Mentions légales du service

Skip to content
Snippets Groups Projects
Commit 5b291966 authored by BESSON Frederic's avatar BESSON Frederic
Browse files

Fix Int63 -> Uint63

parent 2f88542c
No related branches found
Tags 8.13+no
No related merge requests found
...@@ -3,7 +3,7 @@ maintainer: "frederic.besson@inria.fr" ...@@ -3,7 +3,7 @@ maintainer: "frederic.besson@inria.fr"
homepage: "https://gitlab.inria.fr/fbesson/itauto" homepage: "https://gitlab.inria.fr/fbesson/itauto"
dev-repo: "git+https://gitlab.inria.fr/fbesson/itauto.git" dev-repo: "git+https://gitlab.inria.fr/fbesson/itauto.git"
authors: ["Frédéric Besson"] authors: ["Frédéric Besson"]
bug-reports: "frederic.besson@inria.fr" bug-reports: ["frederic.besson@inria.fr" "https://gitlab.inria.fr/fbesson/itauto/-/issues"]
license: "MIT" license: "MIT"
synopsis: "Reflexive SAT solver with Nelson-Oppen support, parameterised by a leaf tactic inside Coq" synopsis: "Reflexive SAT solver with Nelson-Oppen support, parameterised by a leaf tactic inside Coq"
description: """ description: """
...@@ -15,12 +15,16 @@ itauto also provides an SMT-like tactic for propositional reasoning modulo the s ...@@ -15,12 +15,16 @@ itauto also provides an SMT-like tactic for propositional reasoning modulo the s
both arithmetic and function symbols. both arithmetic and function symbols.
""" """
build: [make "-j%{jobs}%"] build: [
[make "-j%{jobs}%"]
[make "test"] {with-test}
]
install: [make "install"] install: [make "install"]
depends: [ depends: [
"ocaml" {>= "4.9~"} "ocaml" {>= "4.9~"}
"coq" {= "dev"} "coq" {= "dev"}
"ocamlbuild" {build} "ocamlbuild" {build}
"coq-mathcomp-zify" {with-test}
] ]
depopts: [ "ocamlformat" {build} ] depopts: [ "ocamlformat" {build} ]
......
...@@ -2,6 +2,7 @@ ...@@ -2,6 +2,7 @@
open Names open Names
open Constr open Constr
module P = ProverPatch module P = ProverPatch
let show_theory_time = let show_theory_time =
......
Require Import Cdcl.Itauto. Require Import Cdcl.Itauto.
Require Import Int63 Bool ZArith Lia. Require Import Uint63 Bool ZArith Lia.
Import Formula. Import Formula.
Import HCons. Import HCons.
......
...@@ -12,7 +12,7 @@ Qed. ...@@ -12,7 +12,7 @@ Qed.
#[local] Instance le_leb : Reflect.RProp2 le := Reflect.mkrProp2 _ _ le leb is_true_le. #[local] Instance le_leb : Reflect.RProp2 le := Reflect.mkrProp2 _ _ le leb is_true_le.
Require Import Cdcl.Itauto. Require Import Cdcl.Itauto.
Require Import Int63. Require Import Uint63.
Lemma map : forall a b, Is_true (a <=? b) -> a <= b. Lemma map : forall a b, Is_true (a <=? b) -> a <= b.
Proof. Proof.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment