2014-08-01 00:48:51 +00:00
|
|
|
----------------------------------------------------------------------------------------------------
|
2014-07-02 14:08:20 +00:00
|
|
|
-- Copyright (c) 2014 Microsoft Corporation. All rights reserved.
|
|
|
|
-- Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
-- Author: Leonardo de Moura
|
2014-08-01 00:48:51 +00:00
|
|
|
----------------------------------------------------------------------------------------------------
|
|
|
|
|
|
|
|
import data.string data.num
|
2014-07-02 02:05:22 +00:00
|
|
|
-- This is just a trick to embed the 'tactic language' as a
|
2014-07-02 14:08:20 +00:00
|
|
|
-- Lean expression. We should view 'tactic' as automation
|
|
|
|
-- that when execute produces a term.
|
2014-09-04 23:36:06 +00:00
|
|
|
-- tactic.builtin is just a "dummy" for creating the
|
2014-07-03 15:06:28 +00:00
|
|
|
-- definitions that are actually implemented in C++
|
2014-07-02 14:08:20 +00:00
|
|
|
inductive tactic : Type :=
|
2014-09-04 23:36:06 +00:00
|
|
|
builtin : tactic
|
|
|
|
|
|
|
|
namespace tactic
|
2014-07-02 02:05:22 +00:00
|
|
|
-- Remark the following names are not arbitrary, the tactic module
|
|
|
|
-- uses them when converting Lean expressions into actual tactic objects.
|
|
|
|
-- The bultin 'by' construct triggers the process of converting a
|
2014-07-02 14:08:20 +00:00
|
|
|
-- a term of type 'tactic' into a tactic that sythesizes a term
|
2014-09-17 21:39:05 +00:00
|
|
|
definition and_then [opaque] (t1 t2 : tactic) : tactic := builtin
|
|
|
|
definition or_else [opaque] (t1 t2 : tactic) : tactic := builtin
|
|
|
|
definition append [opaque] (t1 t2 : tactic) : tactic := builtin
|
|
|
|
definition interleave [opaque] (t1 t2 : tactic) : tactic := builtin
|
|
|
|
definition par [opaque] (t1 t2 : tactic) : tactic := builtin
|
|
|
|
definition fixpoint [opaque] (f : tactic → tactic) : tactic := builtin
|
|
|
|
definition repeat [opaque] (t : tactic) : tactic := builtin
|
|
|
|
definition at_most [opaque] (t : tactic) (k : num) : tactic := builtin
|
|
|
|
definition discard [opaque] (t : tactic) (k : num) : tactic := builtin
|
|
|
|
definition focus_at [opaque] (t : tactic) (i : num) : tactic := builtin
|
|
|
|
definition try_for [opaque] (t : tactic) (ms : num) : tactic := builtin
|
|
|
|
definition now [opaque] : tactic := builtin
|
|
|
|
definition assumption [opaque] : tactic := builtin
|
|
|
|
definition eassumption [opaque] : tactic := builtin
|
|
|
|
definition state [opaque] : tactic := builtin
|
|
|
|
definition fail [opaque] : tactic := builtin
|
|
|
|
definition id [opaque] : tactic := builtin
|
|
|
|
definition beta [opaque] : tactic := builtin
|
|
|
|
definition apply [opaque] {B : Type} (b : B) : tactic := builtin
|
|
|
|
definition unfold [opaque] {B : Type} (b : B) : tactic := builtin
|
|
|
|
definition exact [opaque] {B : Type} (b : B) : tactic := builtin
|
|
|
|
definition trace [opaque] (s : string) : tactic := builtin
|
2014-07-04 17:10:05 +00:00
|
|
|
precedence `;`:200
|
|
|
|
infixl ; := and_then
|
2014-07-03 15:06:28 +00:00
|
|
|
notation `!` t:max := repeat t
|
2014-07-04 17:10:05 +00:00
|
|
|
-- [ t_1 | ... | t_n ] notation
|
|
|
|
notation `[` h:100 `|` r:(foldl 100 `|` (e r, or_else r e) h) `]` := r
|
2014-07-08 21:28:33 +00:00
|
|
|
-- [ t_1 || ... || t_n ] notation
|
|
|
|
notation `[` h:100 `||` r:(foldl 100 `||` (e r, par r e) h) `]` := r
|
2014-07-04 17:10:05 +00:00
|
|
|
definition try (t : tactic) : tactic := [ t | id ]
|
2014-07-03 15:06:28 +00:00
|
|
|
notation `?` t:max := try t
|
2014-07-03 19:59:48 +00:00
|
|
|
definition repeat1 (t : tactic) : tactic := t ; !t
|
|
|
|
definition focus (t : tactic) : tactic := focus_at t 0
|
|
|
|
definition determ (t : tactic) : tactic := at_most t 1
|
2014-08-20 02:32:44 +00:00
|
|
|
|
2014-08-07 23:59:08 +00:00
|
|
|
end tactic
|