Skip to content
GitLab
Projects
Groups
Snippets
/
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in
Toggle navigation
Menu
Open sidebar
Why3
why3
Commits
5619e208
Commit
5619e208
authored
Sep 13, 2015
by
Andrei Paskevich
Browse files
theories/{map,set}.why: remove a warning for map extensionality
parent
ff48ef0d
Changes
2
Hide whitespace changes
Inline
Side-by-side
theories/map.why
View file @
5619e208
...
...
@@ -46,8 +46,10 @@ theory MapExt
predicate (==) (m1 m2: 'a -> 'b) = forall x: 'a. m1 x = m2 x
axiom
extensionality:
lemma
extensionality:
forall m1 m2: 'a -> 'b. m1 == m2 -> m1 = m2
(* This lemma is actually provable in Why3, because of how
eliminate_epsilon handles equality to a lambda-term. *)
end
...
...
theories/set.why
View file @
5619e208
...
...
@@ -129,7 +129,7 @@ theory Set
*)
clone export SetGen with type set = set,
predicate mem = mem,
axiom
extensionality,
predicate mem = mem,
lemma
extensionality,
constant empty = empty, lemma empty_def,
function add = add, lemma add_def,
function remove = remove, lemma remove_def,
...
...
Write
Preview
Supports
Markdown
0%
Try again
or
attach a new file
.
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Cancel
Please
register
or
sign in
to comment