aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-10 14:31:47 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-10 14:31:47 +0000
commitea83ab467124ccdbe2d98434f409a1061b689267 (patch)
tree900d2d2288f5c17184ef80dfb240e841a24dece0 /theories/Structures
parent25533df336888df4255e3882e21d5d5420e5de28 (diff)
Bool: iff lemmas about or, a reflect inductive, an is_true function
For the moment, almost no lemmas about (reflect P b), just the proofs that it is equivalent with an P<->b=true. is_true b is (b=true), and is meant to be added as a coercion if one wants it. In the StdLib, this coercion is not globally activated, but particular files are free to use Local Coercion... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13275 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/Orders.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Structures/Orders.v b/theories/Structures/Orders.v
index d7bdfbf71..f83e77ed8 100644
--- a/theories/Structures/Orders.v
+++ b/theories/Structures/Orders.v
@@ -162,9 +162,9 @@ Module OTF_to_TotalOrder (O:OrderedTypeFull) <: TotalOrder
*)
(** For stating properties like transitivity of [leb],
- we coerce [bool] into [Prop].
- NB: To migrate in Init/Datatype later *)
-Local Coercion is_true b := b = true. (*: bool >-> Sortclass.*)
+ we coerce [bool] into [Prop]. *)
+
+Local Coercion is_true : bool >-> Sortclass.
Hint Unfold is_true.
Module Type HasLeBool (Import T:Typ).