Subject: Ssreflect Users Discussion List
List archive
- From: François Pottier <>
- To:
- Subject: [ssreflect] ssreflect and omega
- Date: Thu, 18 Feb 2016 09:43:17 +0100
Hello,
Once ssreflect is loaded, the tactic "omega" no longer works out of the box
(see attached file for an example). Is there a simple way of expanding away
all of ssreflect's notations and definitions, so that "omega" works again?
Thanks,
--
François Pottier
http://gallium.inria.fr/~fpottier/
Require Import Omega.
Goal
forall x y,
x < y ->
x < y + 1.
Proof.
intros. omega.
Qed.
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq div.
Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
Goal
forall x y,
x < y ->
x < y + 1.
Proof.
intros. omega.
Qed.
- [ssreflect] ssreflect and omega, François Pottier, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Laurent Thery, 02/18/2016
- Re: [ssreflect] ssreflect and omega, François Pottier, 02/18/2016
- Message not available
- Re: [ssreflect] ssreflect and omega, François Pottier, 02/18/2016
- RE: [ssreflect] ssreflect and omega, Georges Gonthier, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Maxime Dénès, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Nicolas Magaud, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Laurent Thery, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Maxime Dénès, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Assia Mahboubi, 02/21/2016
- Re: [ssreflect] ssreflect and omega, François Pottier, 02/22/2016
- Re: [ssreflect] ssreflect and omega, Assia Mahboubi, 02/22/2016
- RE: [ssreflect] ssreflect and omega, Georges Gonthier, 02/18/2016
- Re: [ssreflect] ssreflect and omega, François Pottier, 02/18/2016
- Message not available
- Re: [ssreflect] ssreflect and omega, François Pottier, 02/18/2016
- Re: [ssreflect] ssreflect and omega, Laurent Thery, 02/18/2016
Archive powered by MHonArc 2.6.18.