aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/Depends.thy
blob: d69e663dcc95d90646fbf192982444d7bb9e1e0c (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
(* In order to test the latest thm deps setup, consider this example: *)

theory Depends = Main:

  lemma I: "A ==> A" and K: "A ==> B ==> A" .

(*
This reports I, K depending on several things; for your internal
dependency graph you may interpret this as each member of {I, K} depending
on all the deps.

        Markus
*)

end