aboutsummaryrefslogtreecommitdiff
path: root/lib
diff options
context:
space:
mode:
authorletouzey2010-05-19 15:29:32 +0000
committerletouzey2010-05-19 15:29:32 +0000
commite1feff1215562d8f99fedf73c87011e6d7edca19 (patch)
tree873b23eb1db1430751f3ecb35173d58a0b6a5ff2 /lib
parent6af0706a64f490bea919c39e4a91e09f85c24e23 (diff)
Remove refutpat.ml4, ideal.ml4 is again a normal .ml, let* coded in a naive way
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13017 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'lib')
-rw-r--r--lib/refutpat.ml431
1 files changed, 0 insertions, 31 deletions
diff --git a/lib/refutpat.ml4 b/lib/refutpat.ml4
deleted file mode 100644
index ef28019416..0000000000
--- a/lib/refutpat.ml4
+++ /dev/null
@@ -1,31 +0,0 @@
-(************************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
-(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(************************************************************************)
-
-open Pcaml
-
-(** * Non-irrefutable patterns
-
- This small camlp4 extension creates a "let*" variant of the "let"
- syntax that allow the use of a non-exhaustive pattern. The typical
- usage is:
-
- let* x::l = foo in ...
-
- when foo is already known to be non-empty. This way, no warnings by ocamlc.
- A Failure is raised if the pattern doesn't match the expression.
-*)
-
-
-EXTEND
- expr:
- [[ "let"; "*"; p = patt; "="; e1 = expr; "in"; e2 = expr ->
- <:expr< match $e1$ with
- [ $p$ -> $e2$
- | _ -> failwith "Refutable pattern failed"
- ] >> ]];
-END